src/FOL/ex/.if.thy.ML
author paulson
Thu, 21 Mar 1996 13:02:26 +0100
changeset 1601 0ef6ea27ab15
parent 0 a5a9c433f639
permissions -rw-r--r--
Changes required by removal of the theory argument of Theorem

structure If =
struct

local
 val parse_ast_translation = []
 val parse_preproc = None
 val parse_postproc = None
 val parse_translation = []
 val print_translation = []
 val print_preproc = None
 val print_postproc = None
 val print_ast_translation = []
in

(**** begin of user section ****)

(**** end of user section ****)

val thy = extend_theory (FOL.thy)
 "If"
 ([],
  [],
  [],
  [],
  [(["if"], "[o,o,o]=>o")],
  None)
 [("if_def", "if(P,Q,R) == P&Q | ~P&R")]

val ax = get_axiom thy

val if_def = ax "if_def"


end
end