src/HOL/NumberTheory/Fib.thy
changeset 10147 178deaacb244
parent 9944 2a705d1af4dc
child 11049 7eef34adb852
--- a/src/HOL/NumberTheory/Fib.thy	Tue Oct 03 22:36:22 2000 +0200
+++ b/src/HOL/NumberTheory/Fib.thy	Tue Oct 03 22:37:16 2000 +0200
@@ -6,7 +6,7 @@
 The Fibonacci function.  Demonstrates the use of recdef.
 *)
 
-Fib = Divides + Primes +
+Fib = Primes +
 
 consts fib  :: "nat => nat"
 recdef fib "less_than"