src/HOL/ex/Codegenerator_Pretty.thy
author huffman
Thu, 29 Apr 2010 11:41:04 -0700
changeset 36593 fb69c8cd27bd
parent 31378 d1cbf6393964
permissions -rw-r--r--
define linear algebra concepts using scaleR instead of (op *s); generalized many lemmas, though a few theorems that used to work on type int^'n are a bit less general


(* Author: Florian Haftmann, TU Muenchen *)

header {* Generating code using pretty literals and natural number literals  *}

theory Codegenerator_Pretty
imports "~~/src/HOL/ex/Codegenerator_Candidates" Code_Char Efficient_Nat
begin

declare isnorm.simps [code del]

end