src/HOL/Nominal/Examples/Crary.thy
changeset 22421 51a18dd1ea86
parent 22418 49e2d9744ae1
child 22492 43545e640877
equal deleted inserted replaced
22420:4ccc8c1b08a3 22421:51a18dd1ea86
    29 
    29 
    30 syntax (IfThen output)
    30 syntax (IfThen output)
    31   "==>" :: "prop \<Rightarrow> prop \<Rightarrow> prop"
    31   "==>" :: "prop \<Rightarrow> prop \<Rightarrow> prop"
    32   ("\<^raw:{\rmfamily\upshape\normalsize{}>If\<^raw:\,}> _/ \<^raw:{\rmfamily\upshape\normalsize \,>then\<^raw:\,}>/ _.")
    32   ("\<^raw:{\rmfamily\upshape\normalsize{}>If\<^raw:\,}> _/ \<^raw:{\rmfamily\upshape\normalsize \,>then\<^raw:\,}>/ _.")
    33   "_bigimpl" :: "asms \<Rightarrow> prop \<Rightarrow> prop"
    33   "_bigimpl" :: "asms \<Rightarrow> prop \<Rightarrow> prop"
    34   ("\<^raw:{\rmfamily\upshape\normalsize{}>If\<^raw:\,}> _ /\<^raw:{\rmfamily\upshapce\normalsize \,>then\<^raw:\,}>/ _.")
    34   ("\<^raw:{\rmfamily\upshape\normalsize{}>If\<^raw:\,}> _ /\<^raw:{\rmfamily\upshape\normalsize \,>then\<^raw:\,}>/ _.")
    35   "_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" ("\<^raw:\mbox{>_\<^raw:}> /\<^raw:{\rmfamily\upshape\normalsize \,>and\<^raw:\,}>/ _")
    35   "_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" ("\<^raw:\mbox{>_\<^raw:}> /\<^raw:{\rmfamily\upshape\normalsize \,>and\<^raw:\,}>/ _")
    36   "_asm" :: "prop \<Rightarrow> asms" ("\<^raw:\mbox{>_\<^raw:}>")
    36   "_asm" :: "prop \<Rightarrow> asms" ("\<^raw:\mbox{>_\<^raw:}>")
    37 
    37 
    38 syntax (IfThenNoBox output)
    38 syntax (IfThenNoBox output)
    39   "==>" :: "prop \<Rightarrow> prop \<Rightarrow> prop"
    39   "==>" :: "prop \<Rightarrow> prop \<Rightarrow> prop"