src/HOL/Induct/PropLog.thy
changeset 21404 eb85850d3eb7
parent 20503 503ac4c5ef91
child 23746 a455e69c31cc
--- a/src/HOL/Induct/PropLog.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Induct/PropLog.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -30,7 +30,7 @@
   thms  :: "'a pl set => 'a pl set"
 
 abbreviation
-  thm_rel :: "['a pl set, 'a pl] => bool"   (infixl "|-" 50)
+  thm_rel :: "['a pl set, 'a pl] => bool"   (infixl "|-" 50) where
   "H |- p == p \<in> thms H"
 
 inductive "thms(H)"
@@ -73,7 +73,7 @@
 *}
 
 definition
-  sat :: "['a pl set, 'a pl] => bool"   (infixl "|=" 50)
+  sat :: "['a pl set, 'a pl] => bool"   (infixl "|=" 50) where
     "H |= p  =  (\<forall>tt. (\<forall>q\<in>H. tt[[q]]) --> tt[[p]])"