src/ZF/Induct/PropLog.thy
changeset 24893 b8ef7afe3a6b
parent 20503 503ac4c5ef91
child 35068 544867142ea4
--- a/src/ZF/Induct/PropLog.thy	Sun Oct 07 15:49:25 2007 +0200
+++ b/src/ZF/Induct/PropLog.thy	Sun Oct 07 21:19:31 2007 +0200
@@ -62,8 +62,8 @@
   "is_true_fun(Var(v), t) = (if v \<in> t then 1 else 0)"
   "is_true_fun(p=>q, t) = (if is_true_fun(p,t) = 1 then is_true_fun(q,t) else 1)"
 
-constdefs
-  is_true :: "[i,i] => o"
+definition
+  is_true :: "[i,i] => o"  where
   "is_true(p,t) == is_true_fun(p,t) = 1"
   -- {* this definition is required since predicates can't be recursive *}
 
@@ -84,8 +84,8 @@
   is @{text p}.
 *}
 
-constdefs
-  logcon :: "[i,i] => o"    (infixl "|=" 50)
+definition
+  logcon :: "[i,i] => o"    (infixl "|=" 50)  where
   "H |= p == \<forall>t. (\<forall>q \<in> H. is_true(q,t)) --> is_true(p,t)"