src/HOL/HOL.thy
changeset 17197 917c6e7ca28d
parent 16999 307b2ec590ff
child 17274 746bb4c56800
--- a/src/HOL/HOL.thy	Wed Aug 31 15:46:33 2005 +0200
+++ b/src/HOL/HOL.thy	Wed Aug 31 15:46:34 2005 +0200
@@ -1129,14 +1129,9 @@
   its premise.
 *}
 
-consts
-  "=simp=>" :: "[prop, prop] => prop"  (infixr 1)
-(*
-  "op =simp=>" :: "[prop, prop] => prop"  ("(_/ =simp=> _)" [2, 1] 1)
-syntax
-  "op =simp=>" :: "[prop, prop] => prop"  ("op =simp=>")
-*)
-defs simp_implies_def: "op =simp=> \<equiv> op ==>"
+constdefs
+  simp_implies :: "[prop, prop] => prop"  (infixr "=simp=>" 1)
+  "simp_implies \<equiv> op ==>"
 
 lemma simp_impliesI: 
   assumes PQ: "(PROP P \<Longrightarrow> PROP Q)"